doc-src/Locales/Examples2.thy
changeset 48985 5386df44a037
parent 48984 f51d4a302962
child 48986 037d32448e29
--- a/doc-src/Locales/Examples2.thy	Tue Aug 28 18:46:15 2012 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,24 +0,0 @@
-theory Examples2
-imports Examples
-begin
-text {* \vspace{-5ex} *}
-  interpretation %visible int: partial_order "op \<le> :: [int, int] \<Rightarrow> bool"
-    where "int.less x y = (x < y)"
-  proof -
-    txt {* \normalsize The goals are now:
-      @{subgoals [display]}
-      The proof that~@{text \<le>} is a partial order is as above. *}
-    show "partial_order (op \<le> :: int \<Rightarrow> int \<Rightarrow> bool)"
-      by unfold_locales auto
-    txt {* \normalsize The second goal is shown by unfolding the
-      definition of @{term "partial_order.less"}. *}
-    show "partial_order.less op \<le> x y = (x < y)"
-      unfolding partial_order.less_def [OF `partial_order op \<le>`]
-      by auto
-  qed
-
-text {* Note that the above proof is not in the context of the
-  interpreted locale.  Hence, the premise of @{text
-  "partial_order.less_def"} is discharged manually with @{text OF}.
-  *}
-end