85 lines
3.1 KiB
TeX
85 lines
3.1 KiB
TeX
\documentclass[12pt,a4paper,german]{article}
|
|
\usepackage{url}
|
|
%\usepackage{graphics}
|
|
\usepackage{times}
|
|
\usepackage[T1]{fontenc}
|
|
\usepackage{ngerman}
|
|
\usepackage{float}
|
|
\usepackage{diagbox}
|
|
\usepackage[utf8]{inputenc}
|
|
\usepackage{geometry}
|
|
\usepackage{amsfonts}
|
|
\usepackage{amsmath}
|
|
\usepackage{cancel}
|
|
\usepackage{wasysym}
|
|
\usepackage{csquotes}
|
|
\usepackage{graphicx}
|
|
\usepackage{epsfig}
|
|
\usepackage{paralist}
|
|
\usepackage{tikz}
|
|
\geometry{left=2.0cm,textwidth=17cm,top=3.5cm,textheight=23cm}
|
|
|
|
%%%%%%%%%% Fill out the the definitions %%%%%%%%%
|
|
\def \name {Valentin Brandl} %
|
|
\def \matrikel {108018274494} %
|
|
\def \pname {Marvin Herrmann} %
|
|
\def \pmatrikel {108018265436} %
|
|
\def \gruppe {2 (Mi 10-12 Andre)}
|
|
\def \qname {Pascal Brackmann}
|
|
\def \qmatrikel {108017113834} %
|
|
\def \uebung {7} %
|
|
%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
|
|
|
|
% DO NOT MODIFY THIS HEADER
|
|
\newcommand{\hwsol}{
|
|
\vspace*{-2cm}
|
|
\noindent \matrikel \quad \name \hfill \"Ubungsgruppe: \gruppe \\
|
|
\noindent \pmatrikel \quad \pname \\
|
|
\noindent \qmatrikel \quad \qname \\
|
|
\begin{center}{\Large \bf L\"osung f\"ur \"Ubung \# \uebung}\end{center}
|
|
}
|
|
|
|
\begin{document}
|
|
%Import header
|
|
\hwsol
|
|
|
|
\section*{Aufgabe 7.1}
|
|
|
|
Sei $G=(V,E)$ ein Graph. Mit $G^c := (V,(\frac{V}{2})\setminus E )$ bezeichnen wir den zu G komplementären Graphen. In Hausübung 6.3 wurde definiert, wann ein Graph asymmetrisch ist. Zeige: G ist asymmetrisch $\Leftrightarrow G^c$ ist asymmetrisch\\
|
|
\\
|
|
\noindent
|
|
Definition Asymmetrisch:\\
|
|
Sei $G = (V,E)$ ein ungerichteter Graph. Ein Automorphismus von G ist ein Isomorphismus
|
|
von G auf sich selbst, d.h. eine Bijektion $f : V \rightarrow V$ , so dass $\{u,v\} \in E$ genau dann, wenn
|
|
$\{f(u),f(v)\}g \in E$. Ein Graph heißt genau dann asymmetrisch, wenn die Identität der einzige
|
|
Automorphismus ist.\\
|
|
\\
|
|
\noindent
|
|
\textbf{BEWEIS:}\\
|
|
Seien $G=(V_1,E_1)$ und $G^c=(V_2,E_2)$ zwei Graphen, wobei $G^c$ der Komplementgraph von G ist.\\
|
|
\\
|
|
\noindent
|
|
G hat einen Automorphismus f.\\
|
|
$\Leftrightarrow$\\
|
|
Für alle Kanten $\{u,v\} \in E_1$ ist $\{f(u),f(v)\} \in E_1$ (also eine Kante und gleiches gilt umgekehrt).\\
|
|
$\Leftrightarrow$\\
|
|
Für alle Nichtkanten $\{u,v\} \not \in E_1$ ist $\{f(u),f(v)\} \not \in E_1$ (also keine Kante und gleiches gilt umgekehrt)\\
|
|
$\Leftrightarrow$ (*)(**)\\
|
|
Für alle Kanten $\{u,v\} \in E_2$ ist $\{f(u),f(v)\} \in E_2$ (also eine Kante und gleiches gilt umgekehrt)\\
|
|
$\Leftrightarrow$\\
|
|
Für alle Nichtkanten $\{u,v\} \not \in E_2$ ist $\{f(u),f(v)\} \not \in E_2$ (also keine Kante und gleiches gilt umgekehrt)\\
|
|
$\Leftrightarrow$\\
|
|
$G^c$ hat einen Automorphismus f.\\
|
|
\\
|
|
\noindent
|
|
G asymmetrisch dann ist \textbf{nur} die Identität ein Automorphismus von G und somit auch von $G^c$.
|
|
$G^c$ kann keinen weiteren Automorphismen haben, da dieser sonst einen Automorphismus auf G bildet.\\
|
|
\\
|
|
$G^c$ asymmetrisch dann ist \textbf{nur} die Identität ein Automorphismus von $G^c$ und somit auch von G.
|
|
G kann keinen weiteren Automorphismen haben, da dieser sonst einen Automorphismus auf $G^c$ bildet.\\
|
|
\\
|
|
(*) $\{(u,v)\}$ Kante in G $\Leftrightarrow$ $\{(u,v)\}$ Nichtkante in $G^c$\\
|
|
(**) $\{(u,v)\}$ Nichtkante in G $\Leftrightarrow$ $\{(u,v)\}$ Kante in $G^c$
|
|
|
|
\end{document}
|