src/HOL/HOLCF/Fixrec.thy
changeset 41429 cf5f025bc3c7
parent 41029 f7d8cfa6e7fc
child 42151 4da4fc77664b
equal deleted inserted replaced
41428:44511bf5dcc6 41429:cf5f025bc3c7
   239       (@{const_name spair}, @{const_name match_spair}),
   239       (@{const_name spair}, @{const_name match_spair}),
   240       (@{const_name Pair}, @{const_name match_Pair}),
   240       (@{const_name Pair}, @{const_name match_Pair}),
   241       (@{const_name ONE}, @{const_name match_ONE}),
   241       (@{const_name ONE}, @{const_name match_ONE}),
   242       (@{const_name TT}, @{const_name match_TT}),
   242       (@{const_name TT}, @{const_name match_TT}),
   243       (@{const_name FF}, @{const_name match_FF}),
   243       (@{const_name FF}, @{const_name match_FF}),
   244       (@{const_name UU}, @{const_name match_bottom}) ]
   244       (@{const_name bottom}, @{const_name match_bottom}) ]
   245 *}
   245 *}
   246 
   246 
   247 hide_const (open) succeed fail run
   247 hide_const (open) succeed fail run
   248 
   248 
   249 end
   249 end