Add stuff
All checks were successful
the build was successful

This commit is contained in:
Valentin Brandl 2018-12-04 15:20:35 +01:00
parent c2e3cfa6c7
commit 55f4546a9f
No known key found for this signature in database
GPG Key ID: 30D341DD34118D7D
5 changed files with 96 additions and 26 deletions

View File

@ -0,0 +1,84 @@
\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}

View File

@ -67,10 +67,22 @@
Hamiltonkreis: $(1,3,4,8,10,9,7,5,6,1)$
\begin{figure}[h!]
\centering
\includegraphics[width=0.5\textwidth]{school/di-ma/uebung/07/07_3_b_1.jpg}
\caption{Entfernen eines inneren Knoten}
\end{figure}
\item Entefernen eines äußeren Knoten ($1$):
Hamiltonkreis: $(2,7,9,3,4,5,6,10,8,2)$
\begin{figure}[h!]
\centering
\includegraphics[width=0.5\textwidth]{school/di-ma/uebung/07/07_3_b_2.jpg}
\caption{Entfernen eines äußeren Knoten}
\end{figure}
\end{enumerate}
Für alle (unterscheidbaren) Möglichkeiten, einen Knoten zu entfernen, wurde gezeigt, dass es einen

Binary file not shown.

After

Width:  |  Height:  |  Size: 101 KiB

Binary file not shown.

After

Width:  |  Height:  |  Size: 4.2 MiB

View File

@ -1,26 +0,0 @@
graph {
node [ shape=point ];
1 [ xlabel="1" ];
{
rank="same";
2 [ xlabel="2" ];
}
1 -- 2;
{
rank="same";
3 [ xlabel="3" ];
4 [ xlabel="4" ];
5 [ xlabel="5" ];
6 [ xlabel="6" ];
}
1 -- 3;
1 -- 6;
3 -- 4;
5 -- 6;
7 [ xlabel="7" ];
8 [ xlabel="8" ];
9 [ xlabel="9" ];
10 [ xlabel="10" ];
}