Theory Zippy_Base_Setup

✐‹creator "Kevin Kappelmann"›
chapter ‹Zippy›
theory Zippy_Base_Setup
  imports
    ML_Unification.ML_Logger
    ML_Unification.Setup_Result_Commands
begin

paragraph ‹Summary›
text ‹Zippy is a tree-search framework based on (alternating) zippers.›

setup_result zippy_base_logger = Logger.new_logger Logger.root "Zippy_Base"


end