src/HOL/IOA/meta_theory/Option.ML
changeset 2018 bcd69cc47cf0
parent 2017 dd3e2a91aeca
child 2019 b45d9f2042e0
--- a/src/HOL/IOA/meta_theory/Option.ML	Mon Sep 23 18:26:51 1996 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,23 +0,0 @@
-(*  Title:      Option.ML
-    ID:         $Id$
-    Author:     Tobias Nipkow
-    Copyright   1994  TU Muenchen
-
-Derived rules
-*)
-
-Addsimps [Let_def];
-
-val [prem] = goal Option.thy "P(opt) ==> P(None) | (? x. P(Some(x)))";
- br (prem RS rev_mp) 1;
- by (Option.option.induct_tac "opt" 1);
- by (ALLGOALS(Fast_tac));
-val optE = store_thm("optE", standard(result() RS disjE));
-
-goal Option.thy "x=None | (? y.x=Some(y))"; 
-by (Option.option.induct_tac "x" 1);
-by (Asm_full_simp_tac 1);
-by (rtac disjI2 1);
-by (rtac exI 1);
-by (Asm_full_simp_tac 1);
-qed"opt_cases";