src/HOL/MicroJava/BV/Opt.thy
changeset 12516 d09d0f160888
parent 11085 b830bf10bf71
child 12911 704713ca07ea
--- a/src/HOL/MicroJava/BV/Opt.thy	Sun Dec 16 00:17:18 2001 +0100
+++ b/src/HOL/MicroJava/BV/Opt.thy	Sun Dec 16 00:17:44 2001 +0100
@@ -1,4 +1,4 @@
-(*  Title:      HOL/BCV/Opt.thy
+(*  Title:      HOL/MicroJava/BV/Opt.thy
     ID:         $Id$
     Author:     Tobias Nipkow
     Copyright   2000 TUM
@@ -13,8 +13,8 @@
 constdefs
  le :: "'a ord => 'a option ord"
 "le r o1 o2 == case o2 of None => o1=None |
-                              Some y => (case o1 of None => True |
-                                                    Some x => x <=_r y)"
+                              Some y => (case o1 of None => True
+                                                  | Some x => x <=_r y)"
 
  opt :: "'a set => 'a option set"
 "opt A == insert None {x . ? y:A. x = Some y}"
@@ -22,7 +22,7 @@
  sup :: "'a ebinop => 'a option ebinop"
 "sup f o1 o2 ==  
  case o1 of None => OK o2 | Some x => (case o2 of None => OK o1
-                                              | Some y => (case f x y of Err => Err | OK z => OK (Some z)))"
+     | Some y => (case f x y of Err => Err | OK z => OK (Some z)))"
 
  esl :: "'a esl => 'a option esl"
 "esl == %(A,r,f). (opt A, le r, sup f)"